src/FOLP/ex/If.thy
author wenzelm
Tue, 04 Jul 2006 19:49:54 +0200
changeset 20003 aac2c0d29751
parent 19796 d86e7b1fc472
child 25991 31b38a39e589
permissions -rw-r--r--
polymorphic: always generalize wrt. used_types;

(* $Id$ *)

theory If
imports FOLP
begin

constdefs
  "if" :: "[o,o,o]=>o"
  "if(P,Q,R) == P&Q | ~P&R"

ML {* use_legacy_bindings (the_context ()) *}

end