src/FOLP/ex/If.thy
author wenzelm
Mon, 06 Feb 2006 20:59:11 +0100
changeset 18944 7d2ed9063477
parent 17480 fd19f77dcf60
child 19796 d86e7b1fc472
permissions -rw-r--r--
union_tpairs: Library.merge; Envir.(beta_)eta_contract; tuned;

(* $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