src/FOLP/ex/If.thy
author haftmann
Tue, 10 Jul 2007 17:30:50 +0200
changeset 23709 fd31da8f752a
parent 19796 d86e7b1fc472
child 25991 31b38a39e589
permissions -rw-r--r--
moved lfp_induct2 here
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
17480
fd19f77dcf60 converted to Isar theory format;
wenzelm
parents: 0
diff changeset
     1
(* $Id$ *)
fd19f77dcf60 converted to Isar theory format;
wenzelm
parents: 0
diff changeset
     2
fd19f77dcf60 converted to Isar theory format;
wenzelm
parents: 0
diff changeset
     3
theory If
fd19f77dcf60 converted to Isar theory format;
wenzelm
parents: 0
diff changeset
     4
imports FOLP
fd19f77dcf60 converted to Isar theory format;
wenzelm
parents: 0
diff changeset
     5
begin
fd19f77dcf60 converted to Isar theory format;
wenzelm
parents: 0
diff changeset
     6
fd19f77dcf60 converted to Isar theory format;
wenzelm
parents: 0
diff changeset
     7
constdefs
19796
d86e7b1fc472 quoted "if";
wenzelm
parents: 17480
diff changeset
     8
  "if" :: "[o,o,o]=>o"
17480
fd19f77dcf60 converted to Isar theory format;
wenzelm
parents: 0
diff changeset
     9
  "if(P,Q,R) == P&Q | ~P&R"
fd19f77dcf60 converted to Isar theory format;
wenzelm
parents: 0
diff changeset
    10
fd19f77dcf60 converted to Isar theory format;
wenzelm
parents: 0
diff changeset
    11
ML {* use_legacy_bindings (the_context ()) *}
fd19f77dcf60 converted to Isar theory format;
wenzelm
parents: 0
diff changeset
    12
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    13
end