author | wenzelm |
Wed, 12 Mar 2025 11:39:00 +0100 | |
changeset 82265 | 4b875a4c83b0 |
parent 80914 | d97fdabd9e2b |
permissions | -rw-r--r-- |
62008 | 1 |
(* Title: HOL/HOLCF/IOA/Pred.thy |
40945 | 2 |
Author: Olaf Müller |
17233 | 3 |
*) |
4559 | 4 |
|
62002 | 5 |
section \<open>Logical Connectives lifted to predicates\<close> |
4559 | 6 |
|
17233 | 7 |
theory Pred |
8 |
imports Main |
|
9 |
begin |
|
10 |
||
36452 | 11 |
default_sort type |
4559 | 12 |
|
62005 | 13 |
type_synonym 'a predicate = "'a \<Rightarrow> bool" |
4559 | 14 |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74101
diff
changeset
|
15 |
definition satisfies :: "'a \<Rightarrow> 'a predicate \<Rightarrow> bool" (\<open>_ \<Turnstile> _\<close> [100, 9] 8) |
62005 | 16 |
where "(s \<Turnstile> P) \<longleftrightarrow> P s" |
4559 | 17 |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74101
diff
changeset
|
18 |
definition valid :: "'a predicate \<Rightarrow> bool" (\<open>\<TTurnstile> _\<close> [9] 8) |
62194 | 19 |
where "(\<TTurnstile> P) \<longleftrightarrow> (\<forall>s. (s \<Turnstile> P))" |
4559 | 20 |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74101
diff
changeset
|
21 |
definition Not :: "'a predicate \<Rightarrow> 'a predicate" (\<open>\<^bold>\<not> _\<close> [40] 40) |
74101 | 22 |
where NOT_def: "Not P s \<longleftrightarrow> \<not> P s" |
4559 | 23 |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74101
diff
changeset
|
24 |
definition AND :: "'a predicate \<Rightarrow> 'a predicate \<Rightarrow> 'a predicate" (infixr \<open>\<^bold>\<and>\<close> 35) |
62005 | 25 |
where "(P \<^bold>\<and> Q) s \<longleftrightarrow> P s \<and> Q s" |
4559 | 26 |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74101
diff
changeset
|
27 |
definition OR :: "'a predicate \<Rightarrow> 'a predicate \<Rightarrow> 'a predicate" (infixr \<open>\<^bold>\<or>\<close> 30) |
62005 | 28 |
where "(P \<^bold>\<or> Q) s \<longleftrightarrow> P s \<or> Q s" |
4559 | 29 |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74101
diff
changeset
|
30 |
definition IMPLIES :: "'a predicate \<Rightarrow> 'a predicate \<Rightarrow> 'a predicate" (infixr \<open>\<^bold>\<longrightarrow>\<close> 25) |
62005 | 31 |
where "(P \<^bold>\<longrightarrow> Q) s \<longleftrightarrow> P s \<longrightarrow> Q s" |
4559 | 32 |
|
7661 | 33 |
end |