src/HOL/SMT_Examples/SMT_Examples.thy
changeset 67226 ec32cdaab97b
parent 66758 9312ce5a938d
child 67399 eab6ce8368fa
equal deleted inserted replaced
67225:cb34f5f49a08 67226:ec32cdaab97b
   378   assumes "x * y \<le> 0" and "\<not> y \<le> 0" and "\<not> x \<le> 0"
   378   assumes "x * y \<le> 0" and "\<not> y \<le> 0" and "\<not> x \<le> 0"
   379   shows False
   379   shows False
   380   using assms by (metis mult_le_0_iff)
   380   using assms by (metis mult_le_0_iff)
   381 
   381 
   382 
   382 
   383 subsection {* Linear arithmetic for natural numbers *}
   383 subsection \<open>Linear arithmetic for natural numbers\<close>
   384 
   384 
   385 declare [[smt_nat_as_int]]
   385 declare [[smt_nat_as_int]]
   386 
   386 
   387 lemma "2 * (x::nat) \<noteq> 1" by smt
   387 lemma "2 * (x::nat) \<noteq> 1" by smt
   388 
   388