Skip to main content
Stack Overflow
  1. About
  2. For Teams
Filter by
Sorted by
Tagged with
0 votes
1 answer
109 views

For a uni project I have to create an implication graph from clauses. For example, from the clause (a or b), I can determine these implication : ¬a -> b ¬b -> a but I really can't find the ...
0 votes
2 answers
79 views

I'm new to CPLEX, and I'm doing a project using CP. I have a multilist A that has 4 arguments : one Operation o, one Surgeon s, one Room r and one Time t A[o,s,r,t] == 1 if and only if the operation ...
1 vote
1 answer
470 views

Say I have the following: Lemma my_lemma : forall a b c, a -> (b -> c) -> d. Proof. intros. Then, above the line, I get: X : a X0 : b -> c Let's say that in my proof, I know I'm ...
0 votes
1 answer
239 views

I have just started reading into propositional calculus/logic, and have realised that a lot of the foundational concepts in this area are similar to those encountered in programming. That is, ...
0 votes
2 answers
392 views

Could someone help me linearize this implication? Being x and y integer variables, the implication is the following x >= 1 --> y = 0 y >= 1 --> x = 0 I would really appreciate some help.
0 votes
1 answer
948 views

I have encountered an example property which works here: property p_a; @(posedge clk) $rose(a) -> $rose(b); endproperty There is no syntax error above. Then I tried to modify to this property ...
1 vote
1 answer
155 views

This question is about a project that I am doing, namely, to code Principia Mathematica in Coq. Principia has derived rules of inference, one of which is Syll: ∀ P Q R : Prop, P→Q, Q→R : P→R I am ...
1 vote
1 answer
59 views

Here is a little test: :- begin_tests(tuturuu). test(foo) :- Expected=[a,b],Got=[a,b,c],verdict(foo,Expected,Got). % helper: transform lists A,B into ordered sets As,Bs setify(A,B,As,Bs) :- % ...
4 votes
1 answer
295 views

I see that many theorems in Isabelle/HOL prefer meta-level implication: ==> instead of --> the object logic level, i.e. higher order logic implication. Isabelle wiki says that roughly ...
Gergely's user avatar
  • 7,685
1 vote
1 answer
79 views

Trying to implement and indicator constraint in Python + Gurobi where the indicator(LHS) is a sum of a binary decision variable. Hi, I've would like to implement following in Python + Gurobi: Y_i_d ...
2 votes
1 answer
820 views

I'm trying to prove the transitivity of -> in Coq's propositions: Theorem implies_trans : forall P Q R : Prop, (P -> Q) -> (Q -> R) -> (P -> R). Proof. I wanted to destruct all ...
7 votes
2 answers
1k views

As noted in another StackOverflow answer that I can't seem to find anymore, this pattern emerges frequently in practical Prolog code: pred(X) :- guard(X), ... pred(X) :- \+ guard(X), ....
-1 votes
1 answer
2k views

I'm practicing logical equivalence and I've come across a question that I'm struggling to answer: Show that (R or P -> R or Q) is equivalent to (not R -> (P -> Q)). I've examined the truth tables of ...
-4 votes
1 answer
1k views

I am new into prolog and I've already done some coding, but I have a task I cannot handle. Could you please tell me how to describe a working predicate, that compares arg1, arg2 and arg3 and returns ...
0 votes
1 answer
111 views

I am wondering if there is any way for me to check if a column has a value, if the value is XXXXX then another column must be in the list of (A,B,C). something like: CREATE TABLE test (a CHAR(60),b ...

15 30 50 per page
1
2

AltStyle によって変換されたページ (->オリジナル) /