src/FOL/ex/NewLocaleTest.thy
changeset 29021 ce100fbc3c8e
parent 29019 8e7d6f959bd7
child 29022 54d3a31ca0f6
--- a/src/FOL/ex/NewLocaleTest.thy	Mon Dec 08 14:22:42 2008 +0100
+++ b/src/FOL/ex/NewLocaleTest.thy	Mon Dec 08 18:44:24 2008 +0100
@@ -121,9 +121,14 @@
     and lnot ("-- _" [60] 60)
   assumes assoc: "(x && y) && z = x && (y && z)"
     and notnot: "-- (-- x) = x"
-  defines "x || y == --(-- x && -- y)"
+  defines lor_def: (* FIXME *) "x || y == --(-- x && -- y)"
+begin
 
-print_locale! logic_def
+lemma "x || y = --(-- x && --y)"
+  by (unfold lor_def) (rule refl)
+
+end
+
 
 text {* Theorem statements *}